Skip to content

Commit

Permalink
Require TypingWf in Quotation.ToTemplate.All
Browse files Browse the repository at this point in the history
  • Loading branch information
JasonGross committed Apr 8, 2023
1 parent 554525b commit d2098c0
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions quotation/theories/ToTemplate/All.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
From MetaCoq.Common Require Import config.
From MetaCoq.Template Require Import Ast Typing.
From MetaCoq.Template Require WfAst (*WfTyping*).
From MetaCoq.Quotation.ToTemplate.Template Require Ast Typing WfAst (*WfTyping*).
From MetaCoq.Template Require WfAst TypingWf.
From MetaCoq.Quotation.ToTemplate.Template Require Ast Typing WfAst TypingWf.

(* without typing derivations *)
Module Raw.
Expand All @@ -14,7 +14,7 @@ Module Raw.
Module WfAst.
Definition quote_wf {Σ t} : @WfAst.wf Σ t -> Ast.term := WfAst.quote_wf.
End WfAst.
(* TODO: do we want anything from WfTyping? Is there anything else missing here? *)
(* TODO: do we want anything from TypingWf? Is there anything else missing here? *)
End Raw.

(* eventually we'll have proofs that the above definitions are well-typed *)

0 comments on commit d2098c0

Please sign in to comment.