src/HOL/Library/Case_Converter.thy
changeset 77811 ae9e6218443d
parent 69605 a96320074298
--- 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 \<open>Eliminating pattern matches\<close>
+
 theory Case_Converter
   imports Main
 begin
 
-subsection \<open>Eliminating pattern matches\<close>
-
 definition missing_pattern_match :: "String.literal \<Rightarrow> (unit \<Rightarrow> 'a) \<Rightarrow> 'a" where
   [code del]: "missing_pattern_match m f = f ()"