tuned whitespace;
authorwenzelm
Sun, 27 Dec 2020 17:53:08 +0100
changeset 73015 2d7060a3ea11
parent 73014 90f4df1970b8
child 73016 8644c1efbda2
tuned whitespace;
src/FOL/FOL.thy
src/FOL/IFOL.thy
--- a/src/FOL/FOL.thy	Sun Dec 27 15:55:42 2020 +0100
+++ b/src/FOL/FOL.thy	Sun Dec 27 17:53:08 2020 +0100
@@ -5,8 +5,8 @@
 section \<open>Classical first-order logic\<close>
 
 theory FOL
-imports IFOL
-keywords "print_claset" "print_induct_rules" :: diag
+  imports IFOL
+  keywords "print_claset" "print_induct_rules" :: diag
 begin
 
 ML_file \<open>~~/src/Provers/classical.ML\<close>
--- a/src/FOL/IFOL.thy	Sun Dec 27 15:55:42 2020 +0100
+++ b/src/FOL/IFOL.thy	Sun Dec 27 17:53:08 2020 +0100
@@ -6,8 +6,7 @@
 
 theory IFOL
   imports Pure
-abbrevs "?<" = "\<exists>\<^sub>\<le>\<^sub>1"
-
+  abbrevs "?<" = "\<exists>\<^sub>\<le>\<^sub>1"
 begin
 
 ML_file \<open>~~/src/Tools/misc_legacy.ML\<close>