Skip to content

Commit

Permalink
Merge pull request #108 from buzden/refactor-ttimp-traversals
Browse files Browse the repository at this point in the history
[ refactor ] Compute recursiveness more purely and effectively
  • Loading branch information
buzden authored Mar 28, 2024
2 parents 9bf8554 + 309d67f commit 3b0f6e9
Show file tree
Hide file tree
Showing 6 changed files with 54 additions and 170 deletions.
4 changes: 2 additions & 2 deletions src/Deriving/DepTyCheck/Gen/Checked.idr
Original file line number Diff line number Diff line change
Expand Up @@ -110,7 +110,7 @@ namespace ClojuringCanonicImpl
Yes prf => Just $ Element extSig prf
No _ => Nothing

DerivatorCore => ClojuringContext m => Elaboration m => CanonicGen m where
DerivatorCore => ClojuringContext m => Elaboration m => NamesInfoInTypes => CanonicGen m where
callGen sig fuel values = do

-- check if we are the first, then we need to start the loop
Expand Down Expand Up @@ -172,7 +172,7 @@ namespace ClojuringCanonicImpl
--- Canonic-dischagring function ---

export
runCanonic : DerivatorCore => SortedMap ExternalGenSignature Name -> (forall m. CanonicGen m => m a) -> Elab (a, List Decl)
runCanonic : DerivatorCore => NamesInfoInTypes => SortedMap ExternalGenSignature Name -> (forall m. CanonicGen m => m a) -> Elab (a, List Decl)
runCanonic exts calc = do
let exts = SortedMap.fromList $ exts.asList <&> \namedSig => (fst $ internalise $ fst namedSig, namedSig)
(x, defs, bodies) <- evalRWST exts (empty, empty, True) calc {s=(SortedMap GenSignature Name, List (GenSignature, Name), _)} {w=(_, _)}
Expand Down
6 changes: 3 additions & 3 deletions src/Deriving/DepTyCheck/Gen/Core.idr
Original file line number Diff line number Diff line change
Expand Up @@ -45,10 +45,10 @@ ConstructorDerivator => DerivatorCore where
canonicConsBody sig (consGenName con) con <&> def (consGenName con)

-- calculate which constructors are recursive and which are not
consRecs <- for sig.targetType.cons $ \con => logBounds "consRec" [sig, con] $ do
consRecs <- logBounds "consRec" [sig] $ pure $ sig.targetType.cons <&> \con => do
let conExprs = map type con.args ++ (getExpr <$> snd (unAppAny con.type))
r <- any (hasNameInsideDeep sig.targetType.name) conExprs
pure (con, toRec r)
let r = any (hasNameInsideDeep sig.targetType.name) conExprs
(con, toRec r)

-- decide how to name a fuel argument on the LHS
let fuelArg = "^fuel_arg^" -- I'm using a name containing chars that cannot be present in the code parsed from the Idris frontend
Expand Down
6 changes: 4 additions & 2 deletions src/Deriving/DepTyCheck/Gen/Core/ConsDerive.idr
Original file line number Diff line number Diff line change
Expand Up @@ -37,6 +37,8 @@ namespace NonObligatoryExts
[LeastEffort] {default False simplificationHack : Bool} -> ConstructorDerivator where
consGenExpr sig con givs fuel = do

let niit : NamesInfoInTypes = %search -- I don't why it won't be found without this

-------------------------------------------------------------
-- Prepare intermediate data and functions using this data --
-------------------------------------------------------------
Expand Down Expand Up @@ -114,7 +116,7 @@ namespace NonObligatoryExts
| No _ => fail "INTERNAL ERROR: error in given params set length computation"

-- Check if called subgenerator can call the current one
mutRec <- hasNameInsideDeep sig.targetType.name $ var subsig.targetType.name
let mutRec = hasNameInsideDeep sig.targetType.name $ var subsig.targetType.name

-- Decide whether to use local (decreasing) or outmost fuel, depending on whether we are in mutual recursion with subgen
let subfuel = if mutRec then fuel else var outmostFuelArg
Expand Down Expand Up @@ -159,7 +161,7 @@ namespace NonObligatoryExts
--------------------------------------------------------------------------------

-- Acquire those variables that appear in non-trivial type expressions, i.e. those which needs to be generated before the left-to-right phase
let preLTR = leftToRightArgsTypeApp >>= \(MkTypeApp _ as) => rights (toList as) >>= toList . allVarNames
let preLTR = leftToRightArgsTypeApp >>= \(MkTypeApp _ as) => rights (toList as) >>= allVarNames
let preLTR = SortedSet.fromList $ mapMaybe (flip lookup conArgIdxs) preLTR

-- Find rightmost arguments among `preLTR`
Expand Down
2 changes: 1 addition & 1 deletion src/Deriving/DepTyCheck/Gen/Derive.idr
Original file line number Diff line number Diff line change
Expand Up @@ -44,7 +44,7 @@ Ord GenSignature where
----------------------

public export
interface Elaboration m => CanonicGen m where
interface Elaboration m => NamesInfoInTypes => CanonicGen m where
callGen : (sig : GenSignature) -> (fuel : TTImp) -> Vect sig.givenParams.size TTImp -> m TTImp

export
Expand Down
1 change: 1 addition & 0 deletions src/Deriving/DepTyCheck/Gen/Entry.idr
Original file line number Diff line number Diff line change
Expand Up @@ -296,6 +296,7 @@ deriveGenExpr signature = do
checkResult@(signature ** externals ** _) <- checkTypeIsGen DerivationTask signature
let externalsSigToName = fromList $ externals.externals <&> \(sig, _) => (sig, nameForGen sig)
let fuelArg = outmostFuelArg
niit <- logBounds "namesInfo" [] $ getNamesInfoInTypes signature.targetType
(callExpr, locals) <- runCanonic externalsSigToName $ callMainDerivedGen signature fuelArg
wrapFuel fuelArg <$> internalGenCallingLambda checkResult (local locals callExpr)

Expand Down
205 changes: 43 additions & 162 deletions src/Deriving/DepTyCheck/Util/Reflection.idr
Original file line number Diff line number Diff line change
@@ -1,6 +1,8 @@
||| `Language.Reflection`-related utilities
module Deriving.DepTyCheck.Util.Reflection

import public Control.Applicative.Const

import public Data.Fin
import public Data.Fuel
import public Data.Nat.Pos
Expand Down Expand Up @@ -394,171 +396,50 @@ nameConformsTo cand origin = do

-- simple syntactic search of a `IVar`, disregarding shadowing or whatever
export
allVarNames : TTImp -> LazyList Name
allVarNames expr = ttimp expr where
mutual
allVarNames' : TTImp -> SortedSet Name
allVarNames' = runConst . mapATTImp' f where
f : TTImp -> Const (SortedSet Name) TTImp -> Const (SortedSet Name) TTImp
f (IVar _ n) = const $ MkConst $ singleton n
f _ = id

-- Same as `allVarNames'`, but returning `List`
export
allVarNames : TTImp -> List Name
allVarNames = SortedSet.toList . allVarNames'

export
record NamesInfoInTypes where
constructor Names
names : SortedMap Name $ SortedSet Name

export
hasNameInsideDeep : NamesInfoInTypes => Name -> TTImp -> Bool
hasNameInsideDeep @{tyi} nm = hasInside empty . allVarNames where

ttimp : TTImp -> LazyList Name
ttimp $ IVar _ n = [n]
ttimp $ IPi _ _ z _ argTy retTy = ttimp argTy ++ ttimp retTy ++ piInfo z
ttimp $ ILam _ _ z _ argTy lamTy = ttimp argTy ++ ttimp lamTy ++ piInfo z
ttimp $ ILet _ _ _ _ nTy nVal sc = ttimp nTy ++ ttimp nVal ++ ttimp sc -- should we check `nTy` here?
ttimp $ ICase _ _ _ ty xs = ttimp ty ++ assert_total (foldMap clause xs)
ttimp $ ILocal _ xs y = assert_total (foldMap decl xs) ++ ttimp y
ttimp $ IUpdate _ xs y = assert_total (foldMap fieldUpdate xs) ++ ttimp y
ttimp $ IApp _ y z = ttimp y ++ ttimp z
ttimp $ INamedApp _ y _ w = ttimp y ++ ttimp w
ttimp $ IAutoApp _ y z = ttimp y ++ ttimp z
ttimp $ IWithApp _ y z = ttimp y ++ ttimp z
ttimp $ ISearch _ _ = []
ttimp $ IAlternative _ y xs = altType y ++ assert_total (foldMap ttimp xs)
ttimp $ IRewrite _ y z = ttimp y ++ ttimp z
ttimp $ IBindHere _ _ z = ttimp z
ttimp $ IBindVar _ _ = []
ttimp $ IAs _ _ _ _ w = ttimp w
ttimp $ IMustUnify _ _ z = ttimp z
ttimp $ IDelayed _ _ z = ttimp z
ttimp $ IDelay _ y = ttimp y
ttimp $ IForce _ y = ttimp y
ttimp $ IQuote _ y = ttimp y
ttimp $ IQuoteName _ _ = []
ttimp $ IQuoteDecl _ xs = assert_total $ foldMap decl xs
ttimp $ IUnquote _ y = ttimp y
ttimp $ IPrimVal _ _ = []
ttimp $ IType _ = []
ttimp $ IHole _ _ = []
ttimp $ Implicit _ _ = []
ttimp $ IWithUnambigNames _ _ y = ttimp y

altType : AltType -> LazyList Name
altType FirstSuccess = []
altType Unique = []
altType (UniqueDefault x) = ttimp x

lncpt : List (Name, Count, PiInfo TTImp, TTImp) -> LazyList Name
lncpt = foldMap (\(_, _, pii, tt) => piInfo pii ++ ttimp tt)

ity : ITy -> LazyList Name
ity $ MkTy _ _ _ ty = ttimp ty

decl : Decl -> LazyList Name
decl $ IClaim _ _ _ _ t = ity t
decl $ IData _ _ _ z = data_ z
decl $ IDef _ _ xs = foldMap clause xs
decl $ IParameters _ xs ys = lncpt xs ++ assert_total (foldMap decl ys)
decl $ IRecord _ _ _ _ $ MkRecord _ _ ps _ _ fs = lncpt ps ++ foldMap (\(MkIField _ _ pii _ tt) => piInfo pii ++ ttimp tt) fs
decl $ INamespace _ _ xs = assert_total $ foldMap decl xs
decl $ ITransform _ _ z w = ttimp z ++ ttimp w
decl $ IRunElabDecl _ y = ttimp y
decl $ ILog _ = []
decl $ IBuiltin _ _ _ = []

data_ : Data -> LazyList Name
data_ $ MkData x n tycon _ datacons = maybe [] ttimp tycon ++ foldMap ity datacons
data_ $ MkLater x n tycon = ttimp tycon

fieldUpdate : IFieldUpdate -> LazyList Name
fieldUpdate $ ISetField _ x = ttimp x
fieldUpdate $ ISetFieldApp _ x = ttimp x

clause : Clause -> LazyList Name
clause $ PatClause _ lhs rhs = ttimp lhs ++ ttimp rhs
clause $ WithClause _ lhs _ wval _ _ xs = ttimp lhs ++ ttimp wval ++ assert_total (foldMap clause xs)
clause $ ImpossibleClause _ lhs = ttimp lhs

piInfo : PiInfo TTImp -> LazyList Name
piInfo ImplicitArg = []
piInfo ExplicitArg = []
piInfo AutoImplicit = []
piInfo (DefImplicit x) = ttimp x
hasInside : (visited : SortedSet Name) -> (toLook : List Name) -> Bool
hasInside visited [] = False
hasInside visited (curr::rest) = if curr == nm then True else do
let new = if contains curr visited then [] else maybe [] SortedSet.toList $ lookup curr tyi.names
-- visited is limited and either growing or `new` is empty, thus `toLook` is strictly less
assert_total $ hasInside (insert curr visited) (new ++ rest)

export
hasNameInsideDeep : Elaboration m => Name -> TTImp -> m Bool
hasNameInsideDeep nm expr = evalStateT .| the (SortedSet Name) empty .| hasInside where

hasInside : forall mm. Elaboration mm => MonadState (SortedSet Name) mm => mm Bool
hasInside = ttimp expr where
mutual

ttimp : TTImp -> mm Bool
ttimp $ IVar _ n = if n == nm then pure True else
if contains n !get then pure False else do
modify $ insert n
Just ty <- catch (getInfo' n)
| Nothing => pure False
let subexprs = (map type ty.args) ++ (ty.cons >>= \con => con.type :: map type con.args)
assert_total $ any ttimp subexprs
ttimp $ IPi _ _ z _ argTy retTy = ttimp argTy || ttimp retTy || piInfo z
ttimp $ ILam _ _ z _ argTy lamTy = ttimp argTy || ttimp lamTy || piInfo z
ttimp $ ILet _ _ _ _ nTy nVal sc = ttimp nTy || ttimp nVal || ttimp sc -- should we check `nTy` here?
ttimp $ ICase _ _ _ ty xs = ttimp ty || assert_total (any clause xs)
ttimp $ ILocal _ xs y = assert_total (any decl xs) || ttimp y
ttimp $ IUpdate _ xs y = assert_total (any fieldUpdate xs) || ttimp y
ttimp $ IApp _ y z = ttimp y || ttimp z
ttimp $ INamedApp _ y _ w = ttimp y || ttimp w
ttimp $ IAutoApp _ y z = ttimp y || ttimp z
ttimp $ IWithApp _ y z = ttimp y || ttimp z
ttimp $ ISearch _ _ = pure False
ttimp $ IAlternative _ y xs = altType y || assert_total (any ttimp xs)
ttimp $ IRewrite _ y z = ttimp y || ttimp z
ttimp $ IBindHere _ _ z = ttimp z
ttimp $ IBindVar _ _ = pure False
ttimp $ IAs _ _ _ _ w = ttimp w
ttimp $ IMustUnify _ _ z = ttimp z
ttimp $ IDelayed _ _ z = ttimp z
ttimp $ IDelay _ y = ttimp y
ttimp $ IForce _ y = ttimp y
ttimp $ IQuote _ y = ttimp y
ttimp $ IQuoteName _ _ = pure False
ttimp $ IQuoteDecl _ xs = assert_total $ any decl xs
ttimp $ IUnquote _ y = ttimp y
ttimp $ IPrimVal _ _ = pure False
ttimp $ IType _ = pure False
ttimp $ IHole _ _ = pure False
ttimp $ Implicit _ _ = pure False
ttimp $ IWithUnambigNames _ _ y = ttimp y

altType : AltType -> mm Bool
altType FirstSuccess = pure False
altType Unique = pure False
altType (UniqueDefault x) = ttimp x

lncpt : List (Name, Count, PiInfo TTImp, TTImp) -> mm Bool
lncpt = any (\(_, _, pii, tt) => piInfo pii || ttimp tt)

ity : ITy -> mm Bool
ity $ MkTy _ _ _ ty = ttimp ty

decl : Decl -> mm Bool
decl $ IClaim _ _ _ _ t = ity t
decl $ IData _ _ _ z = data_ z
decl $ IDef _ _ xs = any clause xs
decl $ IParameters _ xs ys = lncpt xs || assert_total (any decl ys)
decl $ IRecord _ _ _ _ $ MkRecord _ _ ps _ _ fs = lncpt ps || any (\(MkIField _ _ pii _ tt) => piInfo pii || ttimp tt) fs
decl $ INamespace _ _ xs = assert_total $ any decl xs
decl $ ITransform _ _ z w = ttimp z || ttimp w
decl $ IRunElabDecl _ y = ttimp y
decl $ ILog _ = pure False
decl $ IBuiltin _ _ _ = pure False

data_ : Data -> mm Bool
data_ $ MkData x n tycon _ datacons = maybe (pure False) ttimp tycon || any ity datacons
data_ $ MkLater x n tycon = ttimp tycon

fieldUpdate : IFieldUpdate -> mm Bool
fieldUpdate $ ISetField _ x = ttimp x
fieldUpdate $ ISetFieldApp _ x = ttimp x

clause : Clause -> mm Bool
clause $ PatClause _ lhs rhs = ttimp lhs || ttimp rhs
clause $ WithClause _ lhs _ wval _ _ xs = ttimp lhs || ttimp wval || assert_total (any clause xs)
clause $ ImpossibleClause _ lhs = ttimp lhs

piInfo : PiInfo TTImp -> mm Bool
piInfo ImplicitArg = pure False
piInfo ExplicitArg = pure False
piInfo AutoImplicit = pure False
piInfo (DefImplicit x) = ttimp x
getNamesInfoInTypes : Elaboration m => TypeInfo -> m NamesInfoInTypes
getNamesInfoInTypes ty = Names <$> go empty [ty]
where

subexprs : TypeInfo -> List TTImp
subexprs ty = map type ty.args ++ (ty.cons >>= \con => con.type :: map type con.args)

go : SortedMap Name (SortedSet Name) -> List TypeInfo -> m $ SortedMap Name $ SortedSet Name
go tyi [] = pure tyi
go tyi (ti::rest) = do
let subes = concatMap allVarNames' $ subexprs ti
new <- map join $ for (SortedSet.toList subes) $ \n =>
if isNothing $ lookup n tyi
then map toList $ catch $ getInfo' n
else pure []
assert_total $ go (insert ti.name subes tyi) (new ++ rest)

public export
isVar : TTImp -> Bool
Expand Down

0 comments on commit 3b0f6e9

Please sign in to comment.