src/Doc/Implementation/Logic.thy
changeset 74266 612b7e0d6721
parent 74200 17090e27aae9
child 74282 c2ee8d993d6a
--- a/src/Doc/Implementation/Logic.thy	Thu Sep 09 10:40:57 2021 +0200
+++ b/src/Doc/Implementation/Logic.thy	Thu Sep 09 12:33:14 2021 +0200
@@ -585,7 +585,7 @@
   @{define_ML Thm.forall_elim: "cterm -> thm -> thm"} \\
   @{define_ML Thm.implies_intr: "cterm -> thm -> thm"} \\
   @{define_ML Thm.implies_elim: "thm -> thm -> thm"} \\
-  @{define_ML Thm.generalize: "Symtab.set * Symtab.set -> int -> thm -> thm"} \\
+  @{define_ML Thm.generalize: "Names.set * Names.set -> int -> thm -> thm"} \\
   @{define_ML Thm.instantiate: "((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list
   -> thm -> thm"} \\
   @{define_ML Thm.add_axiom: "Proof.context ->