# HG changeset patch # User haftmann # Date 1681214342 0 # Node ID ae9e6218443dda4b7da49e5c842d9fd8254f803d # Parent 1a9decb8bfbcf4151e86a53c96a2f97827d642a4 proper section headings diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Cancellation.thy --- a/src/HOL/Library/Cancellation.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Cancellation.thy Tue Apr 11 11:59:02 2023 +0000 @@ -74,7 +74,7 @@ by (auto dest!: le_Suc_ex add_right_imp_eq simp: ab_semigroup_add_class.add_ac(1)) -subsection \Simproc Set-Up\ +text \Simproc Set-Up\ ML_file \Cancellation/cancel.ML\ ML_file \Cancellation/cancel_data.ML\ diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Case_Converter.thy --- a/src/HOL/Library/Case_Converter.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Case_Converter.thy Tue Apr 11 11:59:02 2023 +0000 @@ -1,12 +1,12 @@ (* Author: Pascal Stoop, ETH Zurich Author: Andreas Lochbihler, Digital Asset *) +section \Eliminating pattern matches\ + theory Case_Converter imports Main begin -subsection \Eliminating pattern matches\ - definition missing_pattern_match :: "String.literal \ (unit \ 'a) \ 'a" where [code del]: "missing_pattern_match m f = f ()" diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Code_Cardinality.thy --- a/src/HOL/Library/Code_Cardinality.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Code_Cardinality.thy Tue Apr 11 11:59:02 2023 +0000 @@ -1,4 +1,4 @@ -subsection \Code setup for sets with cardinality type information\ +section \Code setup for sets with cardinality type information\ theory Code_Cardinality imports Cardinality begin diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Code_Test.thy --- a/src/HOL/Library/Code_Test.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Code_Test.thy Tue Apr 11 11:59:02 2023 +0000 @@ -4,6 +4,8 @@ Test infrastructure for the code generator. *) +section \Test infrastructure for the code generator\ + theory Code_Test imports Main keywords "test_code" :: diag diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Extended_Nonnegative_Real.thy --- a/src/HOL/Library/Extended_Nonnegative_Real.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Extended_Nonnegative_Real.thy Tue Apr 11 11:59:02 2023 +0000 @@ -2,7 +2,7 @@ Author: Johannes Hölzl *) -subsection \The type of non-negative extended real numbers\ +section \The type of non-negative extended real numbers\ theory Extended_Nonnegative_Real imports Extended_Real Indicator_Function diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Finite_Lattice.thy --- a/src/HOL/Library/Finite_Lattice.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Finite_Lattice.thy Tue Apr 11 11:59:02 2023 +0000 @@ -2,10 +2,14 @@ Author: Alessandro Coglio *) +section \Finite Lattices\ + theory Finite_Lattice imports Product_Order begin +subsection \Finite Complete Lattices\ + text \A non-empty finite lattice is a complete lattice. Since types are never empty in Isabelle/HOL, a type of classes \<^class>\finite\ and \<^class>\lattice\ diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Lattice_Constructions.thy --- a/src/HOL/Library/Lattice_Constructions.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Lattice_Constructions.thy Tue Apr 11 11:59:02 2023 +0000 @@ -3,12 +3,12 @@ Copyright 2010 TU Muenchen *) +section \Values extended by a bottom element\ + theory Lattice_Constructions imports Main begin -subsection \Values extended by a bottom element\ - datatype 'a bot = Value 'a | Bot instantiation bot :: (preorder) preorder diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Rounded_Division.thy --- a/src/HOL/Library/Rounded_Division.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Rounded_Division.thy Tue Apr 11 11:59:02 2023 +0000 @@ -1,7 +1,7 @@ (* Author: Florian Haftmann, TU Muenchen *) -subsection \Rounded division: modulus centered towards zero.\ +section \Rounded division: modulus centered towards zero.\ theory Rounded_Division imports Main diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Signed_Division.thy --- a/src/HOL/Library/Signed_Division.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Signed_Division.thy Tue Apr 11 11:59:02 2023 +0000 @@ -1,7 +1,7 @@ (* Author: Stefan Berghofer et al. *) -subsection \Signed division: negative results rounded towards zero rather than minus infinity.\ +section \Signed division: negative results rounded towards zero rather than minus infinity.\ theory Signed_Division imports Main