src/Pure/thm.ML
changeset 79270 90c5aadcc4b2
parent 79263 bf2e724ff57e
child 79273 d1e5f6d1ddca
--- a/src/Pure/thm.ML	Sun Dec 17 15:09:55 2023 +0100
+++ b/src/Pure/thm.ML	Sun Dec 17 21:12:18 2023 +0100
@@ -1668,7 +1668,7 @@
               val thy' = Context.certificate_theory cert' handle ERROR msg =>
                 raise CONTEXT (msg, [], [], [th], Option.map Context.Proof opt_ctxt);
 
-              fun zproof p = ZTerm.norm_proof thy' env p;
+              fun zproof p = ZTerm.norm_proof thy' env [full_prop_of th] p;
               fun proof p = Proofterm.norm_proof_remove_types env p;
             in
               Thm (deriv_rule1 zproof proof der,
@@ -2074,7 +2074,7 @@
         val thy' = Context.certificate_theory cert' handle ERROR msg =>
           raise CONTEXT (msg, [], [], [state], Option.map Context.Proof opt_ctxt);
         val normt = Envir.norm_term env;
-        fun zproof p = ZTerm.assumption_proof thy' env Bs Bi n p;
+        fun zproof p = ZTerm.assumption_proof thy' env Bs Bi n [full_prop_of state] p;
         fun proof p =
           Proofterm.assumption_proof (map normt Bs) (normt Bi) n p
           |> not (Envir.is_empty env) ? Proofterm.norm_proof_remove_types env;
@@ -2117,7 +2117,7 @@
     | n =>
         let
           fun zproof p =
-            ZTerm.assumption_proof (Context.certificate_theory cert) Envir.init Bs Bi (n + 1) p;
+            ZTerm.assumption_proof (Context.certificate_theory cert) Envir.init Bs Bi (n + 1) [] p;
           fun proof p = Proofterm.assumption_proof Bs Bi (n + 1) p;
         in
           Thm (deriv_rule1 zproof proof der,
@@ -2371,7 +2371,8 @@
           union_constraints constraints1 constraints2
           |> insert_constraints_env thy' env;
         fun zproof p q =
-          ZTerm.bicompose_proof thy' env smax flatten Bs As A oldAs n (nlift + 1) p q;
+          ZTerm.bicompose_proof thy' env smax flatten Bs As A oldAs n (nlift + 1)
+            [full_prop_of state, full_prop_of orule] p q;
         fun proof p q =
           Proofterm.bicompose_proof env smax flatten Bs As A oldAs n (nlift + 1) p q;
         val th =